Skip to content

Commit

Permalink
test/bugs/github1758.v: add comment explaining tests
Browse files Browse the repository at this point in the history
  • Loading branch information
jdchristensen committed Sep 18, 2023
1 parent 9b9c6d7 commit 5e52ef8
Showing 1 changed file with 2 additions and 0 deletions.
2 changes: 2 additions & 0 deletions test/bugs/github1758.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,8 @@
From HoTT Require Import Basics.Overture HIT.Interval HIT.Flattening Colimits.GraphQuotient
Spaces.Torus.Torus Cubical.

(* Test that various higher inductive types are defined correctly. If they are defined in the most naive way, two uses of the induction principle that are definitionally equal on the point constructors will be considered definitionally equal, which is inconsistent. There is an idiom that must be used in order to force Coq to regard the supplementary data as being required as well. See, for example, Colimits/GraphQuotient.v for the idiom. *)

Fail Definition test_interval (P : interval -> Type) (a : P zero) (b : P one)
(p p' : seg # a = b) :
interval_ind P a b p = interval_ind P a b p'
Expand Down

0 comments on commit 5e52ef8

Please sign in to comment.