View Deliberate.v
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
From mathcomp Require Import ssreflect. | |
Require Import List Nat Ensembles Image. | |
Import ListNotations. | |
Notation empty := (Empty_set _). | |
Notation single := (Singleton _). | |
Notation union := (Union _). | |
Definition bigcup {T} (X : Ensemble (Ensemble T)) : Ensemble T := |
View powcomlat.v
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
From mathcomp Require Import all_ssreflect. | |
Require Import Bool Nat. | |
Set Implicit Arguments. | |
Unset Strict Implicit. | |
Unset Printing Implicit Defensive. | |
Class lattice := Lattice { | |
base : finType; | |
meet : base -> base -> base; |
View OrderLattice.v
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
From mathcomp Require Import all_ssreflect. | |
Require Import Bool. | |
Set Implicit Arguments. | |
Unset Strict Implicit. | |
Unset Printing Implicit Defensive. | |
Class poSet := PoSet { | |
base : finType; |
View Tarski.v
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
From mathcomp Require Export fintype finset ssrbool ssreflect eqtype. | |
Module Type SIG. | |
Parameter T : finType. | |
Parameter A : {set T}. | |
Parameter F : {set T} -> {set T}. | |
Parameter mono : forall (X Y : {set T}), X \subset Y -> F X \subset F Y. | |
End SIG. |
View ArgumentFrame.v
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
From mathcomp Require Export fintype finset ssrbool ssreflect. | |
Module Type FinTypeSig. | |
Parameter T : finType. | |
End FinTypeSig. | |
Module Type ArgFrame (FTS : FinTypeSig). | |
Import FTS. |
View Fixpoint.v
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Require Import Ensembles. | |
From mathcomp Require Import ssreflect. | |
Arguments Singleton {U}. | |
Arguments Union {U}. | |
Arguments Setminus {U}. | |
Arguments Included {U}. | |
Arguments Couple {U}. | |
Arguments Empty_set {U}. |
View resolution.v
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Require Import List Bool Classical. | |
Import ListNotations. | |
From mathcomp Require Import ssreflect ssrbool. | |
Require Import Ensembles ProofIrrelevance Classical_sets. | |
Definition var := nat. | |
Variable fls tru : var. |
View sequent_cal.v
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Require Import List. | |
Import ListNotations. | |
Variable var : Type. | |
Variable tru fls : var. | |
Inductive prop := | |
| Var : var -> prop | |
| Not : prop -> prop | |
| And : prop -> prop -> prop |
View Arguments.v
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
From mathcomp Require Import all_ssreflect. | |
Variables argument position : finType. | |
Definition A := [set : argument]. | |
Definition X := [set : position]. | |
Definition Rel := rel position. | |
Axiom axiomA : 0 < #|argument|. |
View ACTL.v
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Require Export Classical. | |
Module ACTL. | |
Section Def. | |
Context {state action : Set} {trans : state -> action -> state -> Prop} | |
{tau : action} {tau_eq : forall s s', trans s tau s' <-> s = s'}. |
NewerOlder