Theory Ground_Superposition_Example
theory Ground_Superposition_Example
imports
Typed_Ground_Superposition
First_Order_Clause.Monomorphic_Typing
Monomorphic_Superposition
begin
context monomorphic_superposition_calculus
begin
interpretation ground_example: typed_ground_superposition_calculus where
hole = Hole and compose_context = actxt_compose and
apply_context = apply_ground_context and less⇩t = "(≺⇩t⇩G)" and
select = "λ_. {#}" and term_welltyped = "Ground_Term_Typing.welltyped ℱ"
by unfold_locales auto
end
end