TSTP Solution File: SEU221+3 by Drodi---3.5.1

View Problem - Process Solution

%------------------------------------------------------------------------------
% File     : Drodi---3.5.1
% Problem  : SEU221+3 : TPTP v8.1.2. Released v3.2.0.
% Transfm  : none
% Format   : tptp:raw
% Command  : drodi -learnfrom(drodi.lrn) -timeout(%d) %s

% Computer : n004.cluster.edu
% Model    : x86_64 x86_64
% CPU      : Intel(R) Xeon(R) CPU E5-2620 v4 2.10GHz
% Memory   : 8042.1875MB
% OS       : Linux 3.10.0-693.el7.x86_64
% CPULimit : 300s
% WCLimit  : 300s
% DateTime : Wed May 31 12:36:20 EDT 2023

% Result   : Theorem 0.13s 0.37s
% Output   : CNFRefutation 0.13s
% Verified : 
% SZS Type : Refutation
%            Derivation depth      :   11
%            Number of leaves      :   26
% Syntax   : Number of formulae    :  117 (  17 unt;   0 def)
%            Number of atoms       :  434 (  84 equ)
%            Maximal formula atoms :   19 (   3 avg)
%            Number of connectives :  518 ( 201   ~; 209   |;  71   &)
%                                         (  23 <=>;  14  =>;   0  <=;   0 <~>)
%            Maximal formula depth :   18 (   4 avg)
%            Maximal term depth    :    5 (   1 avg)
%            Number of predicates  :   25 (  23 usr;  18 prp; 0-4 aty)
%            Number of functors    :   15 (  15 usr;   4 con; 0-2 aty)
%            Number of variables   :   78 (;  66   !;  12   ?)

% Comments : 
%------------------------------------------------------------------------------
fof(f5,axiom,
    ! [A] :
      ( ( relation(A)
        & function(A) )
     => ( one_to_one(A)
      <=> ! [B,C] :
            ( ( in(B,relation_dom(A))
              & in(C,relation_dom(A))
              & apply(A,B) = apply(A,C) )
           => B = C ) ) ),
    file('/export/starexec/sandbox/benchmark/theBenchmark.p') ).

fof(f6,axiom,
    ! [A] :
      ( ( relation(A)
        & function(A) )
     => ( relation(function_inverse(A))
        & function(function_inverse(A)) ) ),
    file('/export/starexec/sandbox/benchmark/theBenchmark.p') ).

fof(f20,axiom,
    ? [A] :
      ( relation(A)
      & function(A) ),
    file('/export/starexec/sandbox/benchmark/theBenchmark.p') ).

fof(f24,axiom,
    ? [A] :
      ( relation(A)
      & empty(A)
      & function(A) ),
    file('/export/starexec/sandbox/benchmark/theBenchmark.p') ).

fof(f28,axiom,
    ? [A] :
      ( relation(A)
      & function(A)
      & one_to_one(A) ),
    file('/export/starexec/sandbox/benchmark/theBenchmark.p') ).

fof(f35,axiom,
    ! [A] :
      ( ( relation(A)
        & function(A) )
     => ( one_to_one(A)
       => ! [B] :
            ( ( relation(B)
              & function(B) )
           => ( B = function_inverse(A)
            <=> ( relation_dom(B) = relation_rng(A)
                & ! [C,D] :
                    ( ( ( in(C,relation_rng(A))
                        & D = apply(B,C) )
                     => ( in(D,relation_dom(A))
                        & C = apply(A,D) ) )
                    & ( ( in(D,relation_dom(A))
                        & C = apply(A,D) )
                     => ( in(C,relation_rng(A))
                        & D = apply(B,C) ) ) ) ) ) ) ) ),
    file('/export/starexec/sandbox/benchmark/theBenchmark.p') ).

fof(f36,axiom,
    ! [A,B] :
      ( ( relation(B)
        & function(B) )
     => ( ( one_to_one(B)
          & in(A,relation_rng(B)) )
       => ( A = apply(B,apply(function_inverse(B),A))
          & A = apply(relation_composition(function_inverse(B),B),A) ) ) ),
    file('/export/starexec/sandbox/benchmark/theBenchmark.p') ).

fof(f38,conjecture,
    ! [A] :
      ( ( relation(A)
        & function(A) )
     => ( one_to_one(A)
       => one_to_one(function_inverse(A)) ) ),
    file('/export/starexec/sandbox/benchmark/theBenchmark.p') ).

fof(f39,negated_conjecture,
    ~ ! [A] :
        ( ( relation(A)
          & function(A) )
       => ( one_to_one(A)
         => one_to_one(function_inverse(A)) ) ),
    inference(negated_conjecture,[status(cth)],[f38]) ).

fof(f53,plain,
    ! [A] :
      ( ~ relation(A)
      | ~ function(A)
      | ( one_to_one(A)
      <=> ! [B,C] :
            ( ~ in(B,relation_dom(A))
            | ~ in(C,relation_dom(A))
            | apply(A,B) != apply(A,C)
            | B = C ) ) ),
    inference(pre_NNF_transformation,[status(esa)],[f5]) ).

fof(f54,plain,
    ! [A] :
      ( ~ relation(A)
      | ~ function(A)
      | ( ( ~ one_to_one(A)
          | ! [B,C] :
              ( ~ in(B,relation_dom(A))
              | ~ in(C,relation_dom(A))
              | apply(A,B) != apply(A,C)
              | B = C ) )
        & ( one_to_one(A)
          | ? [B,C] :
              ( in(B,relation_dom(A))
              & in(C,relation_dom(A))
              & apply(A,B) = apply(A,C)
              & B != C ) ) ) ),
    inference(NNF_transformation,[status(esa)],[f53]) ).

fof(f55,plain,
    ! [A] :
      ( ~ relation(A)
      | ~ function(A)
      | ( ( ~ one_to_one(A)
          | ! [B,C] :
              ( ~ in(B,relation_dom(A))
              | ~ in(C,relation_dom(A))
              | apply(A,B) != apply(A,C)
              | B = C ) )
        & ( one_to_one(A)
          | ( in(sk0_0(A),relation_dom(A))
            & in(sk0_1(A),relation_dom(A))
            & apply(A,sk0_0(A)) = apply(A,sk0_1(A))
            & sk0_0(A) != sk0_1(A) ) ) ) ),
    inference(skolemization,[status(esa)],[f54]) ).

fof(f57,plain,
    ! [X0] :
      ( ~ relation(X0)
      | ~ function(X0)
      | one_to_one(X0)
      | in(sk0_0(X0),relation_dom(X0)) ),
    inference(cnf_transformation,[status(esa)],[f55]) ).

fof(f58,plain,
    ! [X0] :
      ( ~ relation(X0)
      | ~ function(X0)
      | one_to_one(X0)
      | in(sk0_1(X0),relation_dom(X0)) ),
    inference(cnf_transformation,[status(esa)],[f55]) ).

fof(f59,plain,
    ! [X0] :
      ( ~ relation(X0)
      | ~ function(X0)
      | one_to_one(X0)
      | apply(X0,sk0_0(X0)) = apply(X0,sk0_1(X0)) ),
    inference(cnf_transformation,[status(esa)],[f55]) ).

fof(f60,plain,
    ! [X0] :
      ( ~ relation(X0)
      | ~ function(X0)
      | one_to_one(X0)
      | sk0_0(X0) != sk0_1(X0) ),
    inference(cnf_transformation,[status(esa)],[f55]) ).

fof(f61,plain,
    ! [A] :
      ( ~ relation(A)
      | ~ function(A)
      | ( relation(function_inverse(A))
        & function(function_inverse(A)) ) ),
    inference(pre_NNF_transformation,[status(esa)],[f6]) ).

fof(f62,plain,
    ! [X0] :
      ( ~ relation(X0)
      | ~ function(X0)
      | relation(function_inverse(X0)) ),
    inference(cnf_transformation,[status(esa)],[f61]) ).

fof(f63,plain,
    ! [X0] :
      ( ~ relation(X0)
      | ~ function(X0)
      | function(function_inverse(X0)) ),
    inference(cnf_transformation,[status(esa)],[f61]) ).

fof(f94,plain,
    ( relation(sk0_3)
    & function(sk0_3) ),
    inference(skolemization,[status(esa)],[f20]) ).

fof(f95,plain,
    relation(sk0_3),
    inference(cnf_transformation,[status(esa)],[f94]) ).

fof(f106,plain,
    ( relation(sk0_7)
    & empty(sk0_7)
    & function(sk0_7) ),
    inference(skolemization,[status(esa)],[f24]) ).

fof(f107,plain,
    relation(sk0_7),
    inference(cnf_transformation,[status(esa)],[f106]) ).

fof(f118,plain,
    ( relation(sk0_11)
    & function(sk0_11)
    & one_to_one(sk0_11) ),
    inference(skolemization,[status(esa)],[f28]) ).

fof(f119,plain,
    relation(sk0_11),
    inference(cnf_transformation,[status(esa)],[f118]) ).

fof(f120,plain,
    function(sk0_11),
    inference(cnf_transformation,[status(esa)],[f118]) ).

fof(f138,plain,
    ! [A] :
      ( ~ relation(A)
      | ~ function(A)
      | ~ one_to_one(A)
      | ! [B] :
          ( ~ relation(B)
          | ~ function(B)
          | ( B = function_inverse(A)
          <=> ( relation_dom(B) = relation_rng(A)
              & ! [C,D] :
                  ( ( ~ in(C,relation_rng(A))
                    | D != apply(B,C)
                    | ( in(D,relation_dom(A))
                      & C = apply(A,D) ) )
                  & ( ~ in(D,relation_dom(A))
                    | C != apply(A,D)
                    | ( in(C,relation_rng(A))
                      & D = apply(B,C) ) ) ) ) ) ) ),
    inference(pre_NNF_transformation,[status(esa)],[f35]) ).

fof(f139,plain,
    ! [A,B,C,D] :
      ( pd0_0(D,C,B,A)
    <=> ( ~ in(C,relation_rng(A))
        | D != apply(B,C)
        | ( in(D,relation_dom(A))
          & C = apply(A,D) ) ) ),
    introduced(predicate_definition,[f138]) ).

fof(f140,plain,
    ! [A] :
      ( ~ relation(A)
      | ~ function(A)
      | ~ one_to_one(A)
      | ! [B] :
          ( ~ relation(B)
          | ~ function(B)
          | ( B = function_inverse(A)
          <=> ( relation_dom(B) = relation_rng(A)
              & ! [C,D] :
                  ( pd0_0(D,C,B,A)
                  & ( ~ in(D,relation_dom(A))
                    | C != apply(A,D)
                    | ( in(C,relation_rng(A))
                      & D = apply(B,C) ) ) ) ) ) ) ),
    inference(formula_renaming,[status(thm)],[f138,f139]) ).

fof(f141,plain,
    ! [A] :
      ( ~ relation(A)
      | ~ function(A)
      | ~ one_to_one(A)
      | ! [B] :
          ( ~ relation(B)
          | ~ function(B)
          | ( ( B != function_inverse(A)
              | ( relation_dom(B) = relation_rng(A)
                & ! [C,D] :
                    ( pd0_0(D,C,B,A)
                    & ( ~ in(D,relation_dom(A))
                      | C != apply(A,D)
                      | ( in(C,relation_rng(A))
                        & D = apply(B,C) ) ) ) ) )
            & ( B = function_inverse(A)
              | relation_dom(B) != relation_rng(A)
              | ? [C,D] :
                  ( ~ pd0_0(D,C,B,A)
                  | ( in(D,relation_dom(A))
                    & C = apply(A,D)
                    & ( ~ in(C,relation_rng(A))
                      | D != apply(B,C) ) ) ) ) ) ) ),
    inference(NNF_transformation,[status(esa)],[f140]) ).

fof(f142,plain,
    ! [A] :
      ( ~ relation(A)
      | ~ function(A)
      | ~ one_to_one(A)
      | ! [B] :
          ( ~ relation(B)
          | ~ function(B)
          | ( ( B != function_inverse(A)
              | ( relation_dom(B) = relation_rng(A)
                & ! [C,D] : pd0_0(D,C,B,A)
                & ! [C,D] :
                    ( ~ in(D,relation_dom(A))
                    | C != apply(A,D)
                    | ( in(C,relation_rng(A))
                      & D = apply(B,C) ) ) ) )
            & ( B = function_inverse(A)
              | relation_dom(B) != relation_rng(A)
              | ? [C,D] : ~ pd0_0(D,C,B,A)
              | ? [C,D] :
                  ( in(D,relation_dom(A))
                  & C = apply(A,D)
                  & ( ~ in(C,relation_rng(A))
                    | D != apply(B,C) ) ) ) ) ) ),
    inference(miniscoping,[status(esa)],[f141]) ).

fof(f143,plain,
    ! [A] :
      ( ~ relation(A)
      | ~ function(A)
      | ~ one_to_one(A)
      | ! [B] :
          ( ~ relation(B)
          | ~ function(B)
          | ( ( B != function_inverse(A)
              | ( relation_dom(B) = relation_rng(A)
                & ! [C,D] : pd0_0(D,C,B,A)
                & ! [C,D] :
                    ( ~ in(D,relation_dom(A))
                    | C != apply(A,D)
                    | ( in(C,relation_rng(A))
                      & D = apply(B,C) ) ) ) )
            & ( B = function_inverse(A)
              | relation_dom(B) != relation_rng(A)
              | ~ pd0_0(sk0_14(B,A),sk0_13(B,A),B,A)
              | ( in(sk0_16(B,A),relation_dom(A))
                & sk0_15(B,A) = apply(A,sk0_16(B,A))
                & ( ~ in(sk0_15(B,A),relation_rng(A))
                  | sk0_16(B,A) != apply(B,sk0_15(B,A)) ) ) ) ) ) ),
    inference(skolemization,[status(esa)],[f142]) ).

fof(f144,plain,
    ! [X0,X1] :
      ( ~ relation(X0)
      | ~ function(X0)
      | ~ one_to_one(X0)
      | ~ relation(X1)
      | ~ function(X1)
      | X1 != function_inverse(X0)
      | relation_dom(X1) = relation_rng(X0) ),
    inference(cnf_transformation,[status(esa)],[f143]) ).

fof(f151,plain,
    ! [A,B] :
      ( ~ relation(B)
      | ~ function(B)
      | ~ one_to_one(B)
      | ~ in(A,relation_rng(B))
      | ( A = apply(B,apply(function_inverse(B),A))
        & A = apply(relation_composition(function_inverse(B),B),A) ) ),
    inference(pre_NNF_transformation,[status(esa)],[f36]) ).

fof(f152,plain,
    ! [B] :
      ( ~ relation(B)
      | ~ function(B)
      | ! [A] :
          ( ~ one_to_one(B)
          | ~ in(A,relation_rng(B))
          | ( A = apply(B,apply(function_inverse(B),A))
            & A = apply(relation_composition(function_inverse(B),B),A) ) ) ),
    inference(miniscoping,[status(esa)],[f151]) ).

fof(f153,plain,
    ! [X0,X1] :
      ( ~ relation(X0)
      | ~ function(X0)
      | ~ one_to_one(X0)
      | ~ in(X1,relation_rng(X0))
      | X1 = apply(X0,apply(function_inverse(X0),X1)) ),
    inference(cnf_transformation,[status(esa)],[f152]) ).

fof(f158,plain,
    ? [A] :
      ( relation(A)
      & function(A)
      & one_to_one(A)
      & ~ one_to_one(function_inverse(A)) ),
    inference(pre_NNF_transformation,[status(esa)],[f39]) ).

fof(f159,plain,
    ( relation(sk0_17)
    & function(sk0_17)
    & one_to_one(sk0_17)
    & ~ one_to_one(function_inverse(sk0_17)) ),
    inference(skolemization,[status(esa)],[f158]) ).

fof(f160,plain,
    relation(sk0_17),
    inference(cnf_transformation,[status(esa)],[f159]) ).

fof(f161,plain,
    function(sk0_17),
    inference(cnf_transformation,[status(esa)],[f159]) ).

fof(f162,plain,
    one_to_one(sk0_17),
    inference(cnf_transformation,[status(esa)],[f159]) ).

fof(f163,plain,
    ~ one_to_one(function_inverse(sk0_17)),
    inference(cnf_transformation,[status(esa)],[f159]) ).

fof(f179,plain,
    ! [X0] :
      ( ~ relation(X0)
      | ~ function(X0)
      | ~ one_to_one(X0)
      | ~ relation(function_inverse(X0))
      | ~ function(function_inverse(X0))
      | relation_dom(function_inverse(X0)) = relation_rng(X0) ),
    inference(destructive_equality_resolution,[status(esa)],[f144]) ).

fof(f187,plain,
    ! [X0] :
      ( ~ relation(X0)
      | ~ function(X0)
      | ~ one_to_one(X0)
      | ~ function(function_inverse(X0))
      | relation_dom(function_inverse(X0)) = relation_rng(X0) ),
    inference(forward_subsumption_resolution,[status(thm)],[f179,f62]) ).

fof(f188,plain,
    ( spl0_0
  <=> relation(sk0_17) ),
    introduced(split_symbol_definition) ).

fof(f190,plain,
    ( ~ relation(sk0_17)
    | spl0_0 ),
    inference(component_clause,[status(thm)],[f188]) ).

fof(f191,plain,
    ( spl0_1
  <=> function(sk0_17) ),
    introduced(split_symbol_definition) ).

fof(f193,plain,
    ( ~ function(sk0_17)
    | spl0_1 ),
    inference(component_clause,[status(thm)],[f191]) ).

fof(f194,plain,
    ( spl0_2
  <=> function(function_inverse(sk0_17)) ),
    introduced(split_symbol_definition) ).

fof(f196,plain,
    ( ~ function(function_inverse(sk0_17))
    | spl0_2 ),
    inference(component_clause,[status(thm)],[f194]) ).

fof(f197,plain,
    ( spl0_3
  <=> relation_dom(function_inverse(sk0_17)) = relation_rng(sk0_17) ),
    introduced(split_symbol_definition) ).

fof(f198,plain,
    ( relation_dom(function_inverse(sk0_17)) = relation_rng(sk0_17)
    | ~ spl0_3 ),
    inference(component_clause,[status(thm)],[f197]) ).

fof(f200,plain,
    ( ~ relation(sk0_17)
    | ~ function(sk0_17)
    | ~ function(function_inverse(sk0_17))
    | relation_dom(function_inverse(sk0_17)) = relation_rng(sk0_17) ),
    inference(resolution,[status(thm)],[f187,f162]) ).

fof(f201,plain,
    ( ~ spl0_0
    | ~ spl0_1
    | ~ spl0_2
    | spl0_3 ),
    inference(split_clause,[status(thm)],[f200,f188,f191,f194,f197]) ).

fof(f215,plain,
    ( ~ relation(sk0_17)
    | ~ function(sk0_17)
    | spl0_2 ),
    inference(resolution,[status(thm)],[f196,f63]) ).

fof(f216,plain,
    ( ~ spl0_0
    | ~ spl0_1
    | spl0_2 ),
    inference(split_clause,[status(thm)],[f215,f188,f191,f194]) ).

fof(f218,plain,
    ( $false
    | spl0_1 ),
    inference(forward_subsumption_resolution,[status(thm)],[f193,f161]) ).

fof(f219,plain,
    spl0_1,
    inference(contradiction_clause,[status(thm)],[f218]) ).

fof(f220,plain,
    ( $false
    | spl0_0 ),
    inference(forward_subsumption_resolution,[status(thm)],[f190,f160]) ).

fof(f221,plain,
    spl0_0,
    inference(contradiction_clause,[status(thm)],[f220]) ).

fof(f222,plain,
    ( spl0_6
  <=> relation(function_inverse(sk0_17)) ),
    introduced(split_symbol_definition) ).

fof(f224,plain,
    ( ~ relation(function_inverse(sk0_17))
    | spl0_6 ),
    inference(component_clause,[status(thm)],[f222]) ).

fof(f225,plain,
    ( spl0_7
  <=> one_to_one(function_inverse(sk0_17)) ),
    introduced(split_symbol_definition) ).

fof(f226,plain,
    ( one_to_one(function_inverse(sk0_17))
    | ~ spl0_7 ),
    inference(component_clause,[status(thm)],[f225]) ).

fof(f228,plain,
    ( spl0_8
  <=> in(sk0_1(function_inverse(sk0_17)),relation_rng(sk0_17)) ),
    introduced(split_symbol_definition) ).

fof(f229,plain,
    ( in(sk0_1(function_inverse(sk0_17)),relation_rng(sk0_17))
    | ~ spl0_8 ),
    inference(component_clause,[status(thm)],[f228]) ).

fof(f231,plain,
    ( ~ relation(function_inverse(sk0_17))
    | ~ function(function_inverse(sk0_17))
    | one_to_one(function_inverse(sk0_17))
    | in(sk0_1(function_inverse(sk0_17)),relation_rng(sk0_17))
    | ~ spl0_3 ),
    inference(paramodulation,[status(thm)],[f198,f58]) ).

fof(f232,plain,
    ( ~ spl0_6
    | ~ spl0_2
    | spl0_7
    | spl0_8
    | ~ spl0_3 ),
    inference(split_clause,[status(thm)],[f231,f222,f194,f225,f228,f197]) ).

fof(f233,plain,
    ( spl0_9
  <=> in(sk0_0(function_inverse(sk0_17)),relation_rng(sk0_17)) ),
    introduced(split_symbol_definition) ).

fof(f234,plain,
    ( in(sk0_0(function_inverse(sk0_17)),relation_rng(sk0_17))
    | ~ spl0_9 ),
    inference(component_clause,[status(thm)],[f233]) ).

fof(f236,plain,
    ( ~ relation(function_inverse(sk0_17))
    | ~ function(function_inverse(sk0_17))
    | one_to_one(function_inverse(sk0_17))
    | in(sk0_0(function_inverse(sk0_17)),relation_rng(sk0_17))
    | ~ spl0_3 ),
    inference(paramodulation,[status(thm)],[f198,f57]) ).

fof(f237,plain,
    ( ~ spl0_6
    | ~ spl0_2
    | spl0_7
    | spl0_9
    | ~ spl0_3 ),
    inference(split_clause,[status(thm)],[f236,f222,f194,f225,f233,f197]) ).

fof(f251,plain,
    ( ~ relation(sk0_17)
    | ~ function(sk0_17)
    | spl0_6 ),
    inference(resolution,[status(thm)],[f224,f62]) ).

fof(f252,plain,
    ( ~ spl0_0
    | ~ spl0_1
    | spl0_6 ),
    inference(split_clause,[status(thm)],[f251,f188,f191,f222]) ).

fof(f308,plain,
    ( spl0_23
  <=> one_to_one(sk0_17) ),
    introduced(split_symbol_definition) ).

fof(f310,plain,
    ( ~ one_to_one(sk0_17)
    | spl0_23 ),
    inference(component_clause,[status(thm)],[f308]) ).

fof(f311,plain,
    ( spl0_24
  <=> sk0_1(function_inverse(sk0_17)) = apply(sk0_17,apply(function_inverse(sk0_17),sk0_1(function_inverse(sk0_17)))) ),
    introduced(split_symbol_definition) ).

fof(f312,plain,
    ( sk0_1(function_inverse(sk0_17)) = apply(sk0_17,apply(function_inverse(sk0_17),sk0_1(function_inverse(sk0_17))))
    | ~ spl0_24 ),
    inference(component_clause,[status(thm)],[f311]) ).

fof(f314,plain,
    ( ~ relation(sk0_17)
    | ~ function(sk0_17)
    | ~ one_to_one(sk0_17)
    | sk0_1(function_inverse(sk0_17)) = apply(sk0_17,apply(function_inverse(sk0_17),sk0_1(function_inverse(sk0_17))))
    | ~ spl0_8 ),
    inference(resolution,[status(thm)],[f229,f153]) ).

fof(f315,plain,
    ( ~ spl0_0
    | ~ spl0_1
    | ~ spl0_23
    | spl0_24
    | ~ spl0_8 ),
    inference(split_clause,[status(thm)],[f314,f188,f191,f308,f311,f228]) ).

fof(f317,plain,
    ( $false
    | spl0_23 ),
    inference(forward_subsumption_resolution,[status(thm)],[f310,f162]) ).

fof(f318,plain,
    spl0_23,
    inference(contradiction_clause,[status(thm)],[f317]) ).

fof(f319,plain,
    ( $false
    | ~ spl0_7 ),
    inference(forward_subsumption_resolution,[status(thm)],[f226,f163]) ).

fof(f320,plain,
    ~ spl0_7,
    inference(contradiction_clause,[status(thm)],[f319]) ).

fof(f321,plain,
    ( spl0_25
  <=> sk0_0(function_inverse(sk0_17)) = apply(sk0_17,apply(function_inverse(sk0_17),sk0_0(function_inverse(sk0_17)))) ),
    introduced(split_symbol_definition) ).

fof(f322,plain,
    ( sk0_0(function_inverse(sk0_17)) = apply(sk0_17,apply(function_inverse(sk0_17),sk0_0(function_inverse(sk0_17))))
    | ~ spl0_25 ),
    inference(component_clause,[status(thm)],[f321]) ).

fof(f324,plain,
    ( ~ relation(sk0_17)
    | ~ function(sk0_17)
    | ~ one_to_one(sk0_17)
    | sk0_0(function_inverse(sk0_17)) = apply(sk0_17,apply(function_inverse(sk0_17),sk0_0(function_inverse(sk0_17))))
    | ~ spl0_9 ),
    inference(resolution,[status(thm)],[f234,f153]) ).

fof(f325,plain,
    ( ~ spl0_0
    | ~ spl0_1
    | ~ spl0_23
    | spl0_25
    | ~ spl0_9 ),
    inference(split_clause,[status(thm)],[f324,f188,f191,f308,f321,f233]) ).

fof(f424,plain,
    ( spl0_43
  <=> relation(sk0_11) ),
    introduced(split_symbol_definition) ).

fof(f426,plain,
    ( ~ relation(sk0_11)
    | spl0_43 ),
    inference(component_clause,[status(thm)],[f424]) ).

fof(f427,plain,
    ( spl0_44
  <=> function(sk0_11) ),
    introduced(split_symbol_definition) ).

fof(f429,plain,
    ( ~ function(sk0_11)
    | spl0_44 ),
    inference(component_clause,[status(thm)],[f427]) ).

fof(f443,plain,
    ( spl0_48
  <=> apply(function_inverse(sk0_17),sk0_0(function_inverse(sk0_17))) = apply(function_inverse(sk0_17),sk0_1(function_inverse(sk0_17))) ),
    introduced(split_symbol_definition) ).

fof(f444,plain,
    ( apply(function_inverse(sk0_17),sk0_0(function_inverse(sk0_17))) = apply(function_inverse(sk0_17),sk0_1(function_inverse(sk0_17)))
    | ~ spl0_48 ),
    inference(component_clause,[status(thm)],[f443]) ).

fof(f446,plain,
    ( ~ relation(function_inverse(sk0_17))
    | ~ function(function_inverse(sk0_17))
    | apply(function_inverse(sk0_17),sk0_0(function_inverse(sk0_17))) = apply(function_inverse(sk0_17),sk0_1(function_inverse(sk0_17))) ),
    inference(resolution,[status(thm)],[f59,f163]) ).

fof(f447,plain,
    ( ~ spl0_6
    | ~ spl0_2
    | spl0_48 ),
    inference(split_clause,[status(thm)],[f446,f222,f194,f443]) ).

fof(f461,plain,
    ( spl0_51
  <=> relation(sk0_7) ),
    introduced(split_symbol_definition) ).

fof(f463,plain,
    ( ~ relation(sk0_7)
    | spl0_51 ),
    inference(component_clause,[status(thm)],[f461]) ).

fof(f469,plain,
    ( spl0_53
  <=> relation(sk0_3) ),
    introduced(split_symbol_definition) ).

fof(f471,plain,
    ( ~ relation(sk0_3)
    | spl0_53 ),
    inference(component_clause,[status(thm)],[f469]) ).

fof(f518,plain,
    ( $false
    | spl0_53 ),
    inference(forward_subsumption_resolution,[status(thm)],[f471,f95]) ).

fof(f519,plain,
    spl0_53,
    inference(contradiction_clause,[status(thm)],[f518]) ).

fof(f520,plain,
    ( $false
    | spl0_51 ),
    inference(forward_subsumption_resolution,[status(thm)],[f463,f107]) ).

fof(f521,plain,
    spl0_51,
    inference(contradiction_clause,[status(thm)],[f520]) ).

fof(f522,plain,
    ( $false
    | spl0_44 ),
    inference(forward_subsumption_resolution,[status(thm)],[f429,f120]) ).

fof(f523,plain,
    spl0_44,
    inference(contradiction_clause,[status(thm)],[f522]) ).

fof(f524,plain,
    ( $false
    | spl0_43 ),
    inference(forward_subsumption_resolution,[status(thm)],[f426,f119]) ).

fof(f525,plain,
    spl0_43,
    inference(contradiction_clause,[status(thm)],[f524]) ).

fof(f1019,plain,
    ( spl0_157
  <=> sk0_0(function_inverse(sk0_17)) = sk0_1(function_inverse(sk0_17)) ),
    introduced(split_symbol_definition) ).

fof(f1021,plain,
    ( sk0_0(function_inverse(sk0_17)) != sk0_1(function_inverse(sk0_17))
    | spl0_157 ),
    inference(component_clause,[status(thm)],[f1019]) ).

fof(f1022,plain,
    ( ~ relation(function_inverse(sk0_17))
    | ~ function(function_inverse(sk0_17))
    | sk0_0(function_inverse(sk0_17)) != sk0_1(function_inverse(sk0_17)) ),
    inference(resolution,[status(thm)],[f60,f163]) ).

fof(f1023,plain,
    ( ~ spl0_6
    | ~ spl0_2
    | ~ spl0_157 ),
    inference(split_clause,[status(thm)],[f1022,f222,f194,f1019]) ).

fof(f1031,plain,
    ( sk0_1(function_inverse(sk0_17)) = apply(sk0_17,apply(function_inverse(sk0_17),sk0_0(function_inverse(sk0_17))))
    | ~ spl0_48
    | ~ spl0_24 ),
    inference(backward_demodulation,[status(thm)],[f444,f312]) ).

fof(f1032,plain,
    ( sk0_1(function_inverse(sk0_17)) = sk0_0(function_inverse(sk0_17))
    | ~ spl0_25
    | ~ spl0_48
    | ~ spl0_24 ),
    inference(forward_demodulation,[status(thm)],[f322,f1031]) ).

fof(f1033,plain,
    ( $false
    | spl0_157
    | ~ spl0_25
    | ~ spl0_48
    | ~ spl0_24 ),
    inference(forward_subsumption_resolution,[status(thm)],[f1032,f1021]) ).

fof(f1034,plain,
    ( spl0_157
    | ~ spl0_25
    | ~ spl0_48
    | ~ spl0_24 ),
    inference(contradiction_clause,[status(thm)],[f1033]) ).

fof(f1035,plain,
    $false,
    inference(sat_refutation,[status(thm)],[f201,f216,f219,f221,f232,f237,f252,f315,f318,f320,f325,f447,f519,f521,f523,f525,f1023,f1034]) ).

%------------------------------------------------------------------------------
%----ORIGINAL SYSTEM OUTPUT
% 0.07/0.12  % Problem  : SEU221+3 : TPTP v8.1.2. Released v3.2.0.
% 0.07/0.13  % Command  : drodi -learnfrom(drodi.lrn) -timeout(%d) %s
% 0.13/0.34  % Computer : n004.cluster.edu
% 0.13/0.34  % Model    : x86_64 x86_64
% 0.13/0.34  % CPU      : Intel(R) Xeon(R) CPU E5-2620 v4 @ 2.10GHz
% 0.13/0.34  % Memory   : 8042.1875MB
% 0.13/0.34  % OS       : Linux 3.10.0-693.el7.x86_64
% 0.13/0.34  % CPULimit : 300
% 0.13/0.34  % WCLimit  : 300
% 0.13/0.34  % DateTime : Tue May 30 09:12:52 EDT 2023
% 0.13/0.35  % CPUTime  : 
% 0.13/0.36  % Drodi V3.5.1
% 0.13/0.37  % Refutation found
% 0.13/0.37  % SZS status Theorem for theBenchmark: Theorem is valid
% 0.13/0.37  % SZS output start CNFRefutation for theBenchmark
% See solution above
% 0.13/0.38  % Elapsed time: 0.033399 seconds
% 0.13/0.38  % CPU time: 0.093709 seconds
% 0.13/0.38  % Memory used: 14.154 MB
%------------------------------------------------------------------------------