Skip to content

Commit

Permalink
Use correct scheme kind for CarriersTermAlgebra_ind
Browse files Browse the repository at this point in the history
Elimination is documented as nonrecursive although incorrectly behaves
like Induction until coq/coq#19017
  • Loading branch information
SkySkimmer authored and Alizter committed May 14, 2024
1 parent 23d4007 commit 5a54a54
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion theories/Algebra/Universal/TermAlgebra.v
Original file line number Diff line number Diff line change
Expand Up @@ -30,7 +30,7 @@ Inductive CarriersTermAlgebra {σ} (C : Carriers σ) : Carriers σ :=
DomOperation (CarriersTermAlgebra C) (σ u) ->
CarriersTermAlgebra C (sort_cod (σ u)).

Scheme CarriersTermAlgebra_ind := Elimination for CarriersTermAlgebra Sort Type.
Scheme CarriersTermAlgebra_ind := Induction for CarriersTermAlgebra Sort Type.
Arguments CarriersTermAlgebra_ind {σ}.

Definition CarriersTermAlgebra_rect {σ} := @CarriersTermAlgebra_ind σ.
Expand Down

0 comments on commit 5a54a54

Please sign in to comment.