mirror of
				https://github.com/nmvdw/HITs-Examples
				synced 2025-11-03 23:23:51 +01:00 
			
		
		
		
	Clean up trailing whitespaces and an unused definition.
This commit is contained in:
		@@ -103,21 +103,6 @@ Section operations.
 | 
				
			|||||||
        split ; apply p.
 | 
					        split ; apply p.
 | 
				
			||||||
  Defined.
 | 
					  Defined.
 | 
				
			||||||
 | 
					
 | 
				
			||||||
  Definition map (A B : Type) (f : A -> B) : FSet A -> FSet B.
 | 
					 | 
				
			||||||
  Proof.
 | 
					 | 
				
			||||||
    hrecursion.
 | 
					 | 
				
			||||||
    - apply ∅.
 | 
					 | 
				
			||||||
    - intro a.
 | 
					 | 
				
			||||||
      apply {|f a|}.
 | 
					 | 
				
			||||||
    - apply (∪).
 | 
					 | 
				
			||||||
    - apply assoc.
 | 
					 | 
				
			||||||
    - apply comm.
 | 
					 | 
				
			||||||
    - apply nl.
 | 
					 | 
				
			||||||
    - apply nr.
 | 
					 | 
				
			||||||
    - intros.
 | 
					 | 
				
			||||||
      apply idem.
 | 
					 | 
				
			||||||
  Defined.
 | 
					 | 
				
			||||||
 | 
					 | 
				
			||||||
  Local Ltac remove_transport
 | 
					  Local Ltac remove_transport
 | 
				
			||||||
    := intros ; apply path_forall ; intro Z ; rewrite transport_arrow
 | 
					    := intros ; apply path_forall ; intro Z ; rewrite transport_arrow
 | 
				
			||||||
       ; rewrite transport_const ; simpl.
 | 
					       ; rewrite transport_const ; simpl.
 | 
				
			||||||
 
 | 
				
			|||||||
		Reference in New Issue
	
	Block a user