Skip to content

Commit

Permalink
Fix About info about squashing
Browse files Browse the repository at this point in the history
The previous version is incorrect (it assumes the order is just Prop <= Type with SProp unrelated)
  • Loading branch information
SkySkimmer committed Jun 24, 2024
1 parent 822f40d commit 9d8cf66
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 3 deletions.
4 changes: 2 additions & 2 deletions test-suite/output/Inductive.out
Original file line number Diff line number Diff line change
Expand Up @@ -50,7 +50,7 @@ sempty is universe polymorphic
sempty@{q | } may only be eliminated to produce values whose type is in sort quality q,
unless instantiated such that the quality SProp
is equal to the instantiation of q,
or to Prop or Type if q is instantiated to Type.
or to constant qualities smaller (SProp <= Prop <= Type) than the instantiation of q.
Expands to: Inductive Inductive.sempty
ssig@{q1 q2 q3 | a b} :
forall A : Type@{q1 | a}, (A -> Type@{q2 | b}) -> Type@{q3 | max(a,b)}
Expand All @@ -60,7 +60,7 @@ ssig is universe polymorphic
ssig@{q1 q2 q3 | a b} may only be eliminated to produce values whose type is in sort quality q3,
unless instantiated such that the qualities q1, q2 and Prop
are equal to the instantiation of q3,
or to Prop or Type if q3 is instantiated to Type.
or to constant qualities smaller (SProp <= Prop <= Type) than the instantiation of q3.
Arguments ssig A%type_scope B%function_scope
Expands to: Inductive Inductive.ssig
BoxP@{q | a} : Type@{q | a} -> Prop
Expand Down
2 changes: 1 addition & 1 deletion vernac/prettyp.ml
Original file line number Diff line number Diff line change
Expand Up @@ -240,7 +240,7 @@ let print_squash env ref udecl = match ref with
| QSort (q,_) ->
let ppq = Termops.pr_evd_qvar sigma q in
str "equal to the instantiation of " ++ ppq ++ pr_comma() ++
str "or to Prop or Type if " ++ ppq ++ str " is instantiated to Type"
str "or to constant qualities smaller (SProp <= Prop <= Type) than the instantiation of " ++ ppq
in
let qs = Sorts.Quality.Set.elements qs in
let quality_s, is_s = match qs with
Expand Down

0 comments on commit 9d8cf66

Please sign in to comment.